theory Timed_Automata imports Main begin chapter ‹Basic Definitions and Semantics› section ‹Time› class time = linordered_ab_group_add + assumes dense: "x < y ⟹ ∃z. x < z ∧ z < y" assumes non_trivial: "∃ x. x ≠ 0" begin lemma non_trivial_neg: "∃ x. x < 0" proof - from non_trivial obtain x where "x ≠ 0" by auto then show ?thesis proof (cases "x < 0", auto, goal_cases) case 1 then have "x > 0" by auto then have "(-x) < 0" by auto then show ?case by blast qed qed end