src/HOL/Orderings.thy
changeset 46689 f559866a7aa2
parent 46631 2c5c003cee35
child 46691 72d81e789106
equal deleted inserted replaced
46675:f4ce220d2799 46689:f559866a7aa2
  1297 begin
  1297 begin
  1298 
  1298 
  1299 definition
  1299 definition
  1300   "\<bottom> = (\<lambda>x. \<bottom>)"
  1300   "\<bottom> = (\<lambda>x. \<bottom>)"
  1301 
  1301 
  1302 lemma bot_apply:
  1302 lemma bot_apply (* CANDIDATE [simp, code] *):
  1303   "\<bottom> x = \<bottom>"
  1303   "\<bottom> x = \<bottom>"
  1304   by (simp add: bot_fun_def)
  1304   by (simp add: bot_fun_def)
  1305 
  1305 
  1306 instance proof
  1306 instance proof
  1307 qed (simp add: le_fun_def bot_apply)
  1307 qed (simp add: le_fun_def bot_apply)
  1313 
  1313 
  1314 definition
  1314 definition
  1315   [no_atp]: "\<top> = (\<lambda>x. \<top>)"
  1315   [no_atp]: "\<top> = (\<lambda>x. \<top>)"
  1316 declare top_fun_def_raw [no_atp]
  1316 declare top_fun_def_raw [no_atp]
  1317 
  1317 
  1318 lemma top_apply:
  1318 lemma top_apply (* CANDIDATE [simp, code] *):
  1319   "\<top> x = \<top>"
  1319   "\<top> x = \<top>"
  1320   by (simp add: top_fun_def)
  1320   by (simp add: top_fun_def)
  1321 
  1321 
  1322 instance proof
  1322 instance proof
  1323 qed (simp add: le_fun_def top_apply)
  1323 qed (simp add: le_fun_def top_apply)