merged
authorChristian Urban <urbanc@in.tum.de>
Mon, 15 Feb 2010 17:02:46 +0100
changeset 1156 a6fc645be6e2
parent 1155 5650924c69ed (current diff)
parent 1154 368ec514aa34 (diff)
child 1160 8c65b39bda95
child 1162 6642df770bc4
merged
--- a/Quot/Examples/LarryInt.thy	Mon Feb 15 17:02:26 2010 +0100
+++ b/Quot/Examples/LarryInt.thy	Mon Feb 15 17:02:46 2010 +0100
@@ -1,7 +1,7 @@
 
 header{*The Integers as Equivalence Classes over Pairs of Natural Numbers*}
 
-theory LarryInt 
+theory LarryInt
 imports Nat "../Quotient" "../Quotient_Product"
 begin
 
@@ -373,12 +373,14 @@
   "nat_raw"
 
 abbreviation
-  "less_raw x y \<equiv> (le_raw x y \<and> \<not>(x = y))"
+  "less_raw x y \<equiv> (le_raw x y \<and> \<not>(intrel x y))"
 
 lemma nat_le_eq_zle_raw:
   shows "less_raw (0, 0) w \<or> le_raw (0, 0) z \<Longrightarrow> (nat_raw w \<le> nat_raw z) = (le_raw w z)"
-apply(auto)
-sorry
+  apply (cases w)
+  apply (cases z)
+  apply (simp add: nat_raw_def le_raw_def)
+  by auto
 
 lemma [quot_respect]:
   shows "(intrel ===> op =) nat_raw nat_raw"