diff -r a0c7290a4e27 -r 27cdc0a3a763 Attic/Quot/Examples/IntEx.thy --- a/Attic/Quot/Examples/IntEx.thy Wed Apr 21 12:25:52 2010 +0200 +++ b/Attic/Quot/Examples/IntEx.thy Mon Apr 26 10:01:13 2010 +0200 @@ -165,27 +165,6 @@ apply(lifting plus_assoc_pre) done -lemma int_induct_raw: - assumes a: "P (0::nat, 0)" - and b: "\i. P i \ P (my_plus i (1,0))" - and c: "\i. P i \ P (my_plus i (my_neg (1,0)))" - shows "P x" - apply(case_tac x) apply(simp) - apply(rule_tac x="b" in spec) - apply(rule_tac Nat.induct) - apply(rule allI) - apply(rule_tac Nat.induct) - using a b c apply(auto) - done - -lemma int_induct: - assumes a: "P ZERO" - and b: "\i. P i \ P (PLUS i ONE)" - and c: "\i. P i \ P (PLUS i (NEG ONE))" - shows "P x" - using a b c - by (lifting int_induct_raw) - lemma ex1tst: "Bex1_rel (op \) (\x :: nat \ nat. x \ x)" sorry