# HG changeset patch # User huffman # Date 1288219801 25200 # Node ID b5e1ab22198aeb059a381b10c333fa9d15db8caa # Parent 4cce7c7084027360ac2673260f3d92f1459165ea rename constant trifte to tr_case diff -r 4cce7c708402 -r b5e1ab22198a src/HOLCF/Tr.thy --- a/src/HOLCF/Tr.thy Wed Oct 27 14:31:39 2010 -0700 +++ b/src/HOLCF/Tr.thy Wed Oct 27 15:50:01 2010 -0700 @@ -64,24 +64,23 @@ default_sort pcpo -definition - trifte :: "'c \ 'c \ tr \ 'c" where - ifte_def: "trifte = (\ t e. FLIFT b. if b then t else e)" +definition tr_case :: "'a \ 'a \ tr \ 'a" where + "tr_case = (\ t e (Def b). if b then t else e)" abbreviation cifte_syn :: "[tr, 'c, 'c] \ 'c" ("(If (_)/ then (_)/ else (_))" [0, 0, 60] 60) where - "If b then e1 else e2 == trifte\e1\e2\b" + "If b then e1 else e2 == tr_case\e1\e2\b" translations - "\ (XCONST TT). t" == "CONST trifte\t\\" - "\ (XCONST FF). t" == "CONST trifte\\\t" + "\ (XCONST TT). t" == "CONST tr_case\t\\" + "\ (XCONST FF). t" == "CONST tr_case\\\t" lemma ifte_thms [simp]: "If \ then e1 else e2 = \" "If FF then e1 else e2 = e2" "If TT then e1 else e2 = e1" -by (simp_all add: ifte_def TT_def FF_def) +by (simp_all add: tr_case_def TT_def FF_def) subsection {* Boolean connectives *} @@ -110,7 +109,7 @@ text {* tactic for tr-thms with case split *} -lemmas tr_defs = andalso_def orelse_def neg_def ifte_def TT_def FF_def +lemmas tr_defs = andalso_def orelse_def neg_def tr_case_def TT_def FF_def text {* lemmas about andalso, orelse, neg and if *}