changeset 195 | 72165b83b9d6 |
parent 194 | 03c03e88efa9 |
parent 193 | b888119a18ff |
child 196 | 9163c0f9830d |
--- a/IntEx.thy Mon Oct 26 15:31:53 2009 +0100 +++ b/IntEx.thy Mon Oct 26 15:32:17 2009 +0100 @@ -23,6 +23,13 @@ term ZERO thm ZERO_def +(* +quotient_def (with my_int) + ZERO :: "my_int" +where + "ZERO \<equiv> (0::nat, 0::nat)" +*) + local_setup {* make_const_def @{binding ONE} @{term "(1::nat, 0::nat)"} NoSyn @{typ "nat \<times> nat"} @{typ "my_int"} #> snd *}